src/HOL/Bali/DefiniteAssignment.thy
changeset 72610 00fce84413db
parent 69597 ff784d5a5bfb
child 77645 7edbb16bc60f
--- a/src/HOL/Bali/DefiniteAssignment.thy	Sun Nov 15 13:06:41 2020 +0000
+++ b/src/HOL/Bali/DefiniteAssignment.thy	Sun Nov 15 13:08:13 2020 +0000
@@ -566,7 +566,7 @@
      in this rule. For example, if \<^term>\<open>e\<close> is constantly \<^term>\<open>True\<close> then 
      \<^term>\<open>assigns_if False e = UNIV\<close> and therefor \<^term>\<open>nrm C2=UNIV\<close>.
      So finally \<^term>\<open>nrm A = nrm C1\<close>. For the break maps this trick 
-     workd too, because the trival break map will map all labels to 
+     workd too, because the trivial break map will map all labels to 
      \<^term>\<open>UNIV\<close>. In the example, if no break occurs in \<^term>\<open>c2\<close> the break
      maps will trivially map to \<^term>\<open>UNIV\<close> and if a break occurs it will map
      to \<^term>\<open>UNIV\<close> too, because \<^term>\<open>assigns_if False e = UNIV\<close>. So