Admin/polyml/future/run
author bulwahn
Tue, 08 May 2012 14:31:03 +0200
changeset 47893 4cf901b1089a
parent 44155 ae2906662eec
permissions -rwxr-xr-x
specialised fact in the Record theory should not be appear in proofs discovered by sledgehammer
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
44153
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     1
#!/bin/bash
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     2
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     3
POLY="${1:-poly}"
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     4
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     5
THIS="$(cd $(dirname "$0"); pwd)"
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     6
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     7
cd "$THIS/../../../src/Pure"
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
     8
echo "use \"../../Admin/polyml/future/ROOT.ML\";"
44155
wenzelm
parents: 44153
diff changeset
     9
exec "$POLY"
44153
aefbb5cc8908 minimal script to run raw Poly/ML with concurrency library;
wenzelm
parents:
diff changeset
    10