- Set your
XCURSOR_SIZE
to 32 (or desired size) in either your/etc/nixos/configuration.nix
environment.variables.XCURSOR_SIZE = "32";
or ~/.Xresources
:
@Iceland_jack: https://twitter.com/Iceland_jack/status/1130243968820830208 | |
< begin :: ([a] -> res) -> res | |
< begin k = k [] | |
< push :: [a] -> a -> ([a] -> res) -> res | |
< push as a k = k (a : as) | |
< add :: Num a => [a] -> ([a] -> res) -> res | |
< add (a:b:rest) k = k (b+a:rest) |
{-# LANGUAGE DeriveFunctor #-} | |
import Control.Arrow ((&&&)) | |
import Data.Bifunctor | |
-- Recursion Schemes for Dynamic Programming | |
-- Kabanov and Vene, Mathematics for Program Construction 2006 | |
-- Basic stuff | |
newtype Mu f = In { out :: f (Mu f) } |
{-# LANGUAGE ExistentialQuantification, RankNTypes #-} | |
module Main where | |
{-@ LIQUID "--higherorder" @-} | |
import Language.Haskell.Liquid.ProofCombinators | |
import Data.Functor.Const | |
import Data.Functor.Identity | |
type Lens s t a b = forall f. Functor f => (a -> f b) -> (s -> f t) |
{-# LANGUAGE | |
DataKinds | |
, TypeApplications | |
, TypeFamilies | |
, TypeOperators | |
, TypeInType | |
, KindSignatures | |
, ExistentialQuantification | |
, InstanceSigs | |
, ScopedTypeVariables |
Require Import Coq.Lists.List. | |
Open Scope bool_scope. | |
(* This is a direct definition of CGTs, using just one inductive type | |
instead of a pair of mutually-inductive types *) | |
Inductive game := Game { | |
left_moves : list game; | |
right_moves : list game |
{-# LANGUAGE FlexibleInstances #-} | |
-- | Fun with typeclasses | |
module Box where | |
import Prelude hiding (Functor(..), Applicative(..), Monad(..), Monoid(..), (.)) | |
infixr 6 <> | |
-------------------------------------------------------------------------------- | |
-- * Parametricity and typeclasses | |
-- see https://www.schoolofhaskell.com/school/starting-with-haskell/introduction-to-haskell/5-type-classes |
gnuindent -kr -l80 -ut -i8 -ts8 -sob *.c *.h | |
# cribbed from scripts/Lindent from kernel | |
gnuindent -npro -kr -i8 -ts8 -sob -l80 -ss -ncs -cp1 |
#! /usr/bin/runhaskell | |
{-# LANGUAGE FlexibleContexts #-} | |
module Lib where | |
import Diagrams.Prelude | |
import Diagrams.Backend.PGF.CmdLine | |
pipeline :: Diagram PGF | |
pipeline = foldr1 (|||) labelledBlocks | |
where |
I hereby claim:
To claim this, I am signing this object: