src/HOL/HOL.thy
changeset 41229 d797baa3d57c
parent 41184 5c6f44d22f51
child 41251 1e6d86821718
--- a/src/HOL/HOL.thy	Fri Dec 17 17:08:56 2010 +0100
+++ b/src/HOL/HOL.thy	Fri Dec 17 17:43:54 2010 +0100
@@ -103,9 +103,8 @@
 notation (xsymbols)
   iff  (infixr "\<longleftrightarrow>" 25)
 
-nonterminals
-  letbinds  letbind
-  case_syn  cases_syn
+nonterminal letbinds and letbind
+nonterminal case_syn and cases_syn
 
 syntax
   "_The"        :: "[pttrn, bool] => 'a"                 ("(3THE _./ _)" [0, 10] 10)