src/HOL/HOL.thy
changeset 41251 1e6d86821718
parent 41247 c5cb19ecbd41
parent 41229 d797baa3d57c
child 41636 934b4ad9b611
equal deleted inserted replaced
41247:c5cb19ecbd41 41251:1e6d86821718
   101   "A <-> B == A = B"
   101   "A <-> B == A = B"
   102 
   102 
   103 notation (xsymbols)
   103 notation (xsymbols)
   104   iff  (infixr "\<longleftrightarrow>" 25)
   104   iff  (infixr "\<longleftrightarrow>" 25)
   105 
   105 
   106 nonterminals
   106 nonterminal letbinds and letbind
   107   letbinds  letbind
   107 nonterminal case_syn and cases_syn
   108   case_syn  cases_syn
       
   109 
   108 
   110 syntax
   109 syntax
   111   "_The"        :: "[pttrn, bool] => 'a"                 ("(3THE _./ _)" [0, 10] 10)
   110   "_The"        :: "[pttrn, bool] => 'a"                 ("(3THE _./ _)" [0, 10] 10)
   112 
   111 
   113   "_bind"       :: "[pttrn, 'a] => letbind"              ("(2_ =/ _)" 10)
   112   "_bind"       :: "[pttrn, 'a] => letbind"              ("(2_ =/ _)" 10)