src/HOL/HOL.thy
changeset 62521 6383440f41a8
parent 62390 842917225d56
child 62522 d32c23d29968
equal deleted inserted replaced
62520:2382876c238b 62521:6383440f41a8
   153 notation (ASCII)
   153 notation (ASCII)
   154   All  (binder "ALL " 10) and
   154   All  (binder "ALL " 10) and
   155   Ex  (binder "EX " 10) and
   155   Ex  (binder "EX " 10) and
   156   Ex1  (binder "EX! " 10)
   156   Ex1  (binder "EX! " 10)
   157 
   157 
   158 notation (HOL)
   158 notation (input)
   159   All  (binder "! " 10) and
   159   All  (binder "! " 10) and
   160   Ex  (binder "? " 10) and
   160   Ex  (binder "? " 10) and
   161   Ex1  (binder "?! " 10)
   161   Ex1  (binder "?! " 10)
   162 
   162 
   163 
   163