File tree 3 files changed +4
-2
lines changed
3 files changed +4
-2
lines changed Original file line number Diff line number Diff line change @@ -134,8 +134,10 @@ sizedTypesModules = map modToFile
134
134
, " Data.Container.Any"
135
135
, " Data.Container.FreeMonad"
136
136
, " Data.Nat.PseudoRandom.LCG.Unsafe"
137
+ , " Data.Tree.Binary.Show"
137
138
, " Data.Tree.Rose"
138
139
, " Data.Tree.Rose.Properties"
140
+ , " Data.Tree.Rose.Show"
139
141
, " Data.Trie"
140
142
, " Data.Trie.NonEmpty"
141
143
, " Relation.Unary.Sized"
Original file line number Diff line number Diff line change 4
4
-- 1 dimensional pretty printing of binary trees
5
5
------------------------------------------------------------------------
6
6
7
- {-# OPTIONS --without-K --safe -- sized-types #-}
7
+ {-# OPTIONS --without-K --sized-types #-}
8
8
9
9
open import Level using (Level)
10
10
open import Data.List.Base as List using (List; []; [_]; _∷_; _∷ʳ_)
Original file line number Diff line number Diff line change 4
4
-- 1 dimensional pretty printing of rose trees
5
5
------------------------------------------------------------------------
6
6
7
- {-# OPTIONS --without-K --safe -- sized-types #-}
7
+ {-# OPTIONS --without-K --sized-types #-}
8
8
9
9
module Data.Tree.Rose.Show where
10
10
You can’t perform that action at this time.
0 commit comments